Skip to content

Commit

Permalink
use inline ring solver
Browse files Browse the repository at this point in the history
  • Loading branch information
mzeuner committed Feb 26, 2024
1 parent 9f02434 commit e582d07
Showing 1 changed file with 1 addition and 4 deletions.
5 changes: 1 addition & 4 deletions Cubical/Algebra/ZariskiLattice/Properties.agda
Original file line number Diff line number Diff line change
Expand Up @@ -101,11 +101,8 @@ module _ (R : CommRing ℓ) where
f ∈ₚ R ˣ
fgHelper (α , 1ⁿ≡α₀f+0) = α zero , path
where
useSolver : f α₀ f · α₀ ≡ α₀ · f + 0r
useSolver = solve R

path : f · α zero ≡ 1r
path = f · α zero ≡⟨ useSolver _ _
path = f · α zero ≡⟨ solve! R
α zero · f + 0r ≡⟨ sym 1ⁿ≡α₀f+0 ⟩
1r ^ n ≡⟨ 1ⁿ≡1 n ⟩
1r ∎
Expand Down

0 comments on commit e582d07

Please sign in to comment.