Skip to content

Commit

Permalink
Fix typo
Browse files Browse the repository at this point in the history
Signed-off-by: Sky Wilshaw <zeramorphic@proton.me>
  • Loading branch information
zeramorphic committed Oct 27, 2024
1 parent 2b3abe8 commit 5c54e26
Showing 1 changed file with 2 additions and 2 deletions.
4 changes: 2 additions & 2 deletions ConNF/Counting/Strong.lean
Original file line number Diff line number Diff line change
Expand Up @@ -180,7 +180,7 @@ def preStrong (S : Support β) : Support β :=

theorem le_preStrong (S : Support β) :
S ≤ S.preStrong :=
le_add.trans le_add
le_add_right.trans le_add_right

theorem preStrong_atoms (S : Support β) (A : β ↝ ⊥) :
(S.preStrong ⇘. A)ᴬ = (S ⇘. A)ᴬ + ((S + S.constrainsNearLitters).constrainsAtoms ⇘. A)ᴬ := by
Expand Down Expand Up @@ -243,7 +243,7 @@ def strong (S : Support β) : Support β :=

theorem preStrong_le_strong (S : Support β) :
S.preStrong ≤ S.strong :=
le_add
le_add_right

theorem le_strong (S : Support β) :
S ≤ S.strong :=
Expand Down

0 comments on commit 5c54e26

Please sign in to comment.