Skip to content

Commit

Permalink
Some updates
Browse files Browse the repository at this point in the history
Signed-off-by: zeramorphic <[email protected]>
  • Loading branch information
zeramorphic committed Oct 24, 2024
1 parent a2b708e commit 122b11a
Show file tree
Hide file tree
Showing 4 changed files with 284 additions and 22 deletions.
4 changes: 4 additions & 0 deletions ConNF/Aux/Rel.lean
Original file line number Diff line number Diff line change
Expand Up @@ -80,6 +80,10 @@ theorem codomEqDom_iff' (r : Rel α α) :
theorem OneOne.inv {r : Rel α β} (h : r.OneOne) : r.inv.OneOne :=
⟨⟨h.coinjective⟩, ⟨h.injective⟩⟩

theorem inv_apply {r : Rel α β} {x : α} {y : β} :
r.inv y x ↔ r x y :=
Iff.rfl

theorem inv_injective : Function.Injective (inv : Rel α β → Rel β α) := by
intro r s h
ext a b : 2
Expand Down
21 changes: 18 additions & 3 deletions ConNF/Counting/CodingFunction.lean
Original file line number Diff line number Diff line change
Expand Up @@ -87,13 +87,13 @@ theorem ext_aux {χ₁ χ₂ : CodingFunction β} {S : Support β} {x : TSet β}
exact χ₂.smul_rel h₂ ρ

theorem ext {χ₁ χ₂ : CodingFunction β} (S : Support β) (x : TSet β)
(h : χ₁.rel S x χ₂.rel S x) :
(h : χ₁.rel S x) (h₂ : χ₂.rel S x) :
χ₁ = χ₂ := by
apply ext'
intro _ _
constructor
· apply ext_aux h.1 h.2
· apply ext_aux h.2 h.1
· apply ext_aux h₁ h₂
· apply ext_aux h₂ h₁

end CodingFunction

Expand Down Expand Up @@ -122,4 +122,19 @@ theorem Tangle.code_rel_self (t : Tangle β) :
use 1
simp only [allPermForget_one, one_smul, and_self]

theorem Tangle.code_eq_code_iff (t₁ t₂ : Tangle β) :
t₁.code = t₂.code ↔ ∃ ρ : AllPerm β, ρ • t₁ = t₂ := by
constructor
· intro h
have := t₂.code_rel_self
rw [← h] at this
obtain ⟨ρ, hρ₁, hρ₂⟩ := this
use ρ
exact Tangle.ext hρ₂ hρ₁
· rintro ⟨ρ, rfl⟩
symm
apply CodingFunction.ext _ _ (ρ • t₁).code_rel_self
use ρ
exact ⟨rfl, rfl⟩

end ConNF
Loading

0 comments on commit 122b11a

Please sign in to comment.