Documentation

ConNF.Model.ConstructHypothesis

New file #

In this file...

Main declarations #

def ConNF.constructAllPermSderiv [Params] {α : Λ} (M : (β : Λ) → β < αMotive β) (H : (β : Λ) → (h : β < α) → Hypothesis (M β h) fun (γ : Λ) (h' : γ < β) => M γ ) {β : Λ} (h : β < α) (ρ : AllPerm α) :
AllPerm β
Equations
Instances For
    def ConNF.constructAllPermBotSderiv [Params] {α : Λ} (M : (β : Λ) → β < αMotive β) (H : (β : Λ) → (h : β < α) → Hypothesis (M β h) fun (γ : Λ) (h' : γ < β) => M γ ) (ρ : AllPerm α) :
    Equations
    Instances For
      def ConNF.constructSingleton [Params] {α : Λ} (M : (β : Λ) → β < αMotive β) (H : (β : Λ) → (h : β < α) → Hypothesis (M β h) fun (γ : Λ) (h' : γ < β) => M γ ) {β : Λ} (h : β < α) (x : TSet β) :
      TSet α
      Equations
      Instances For
        theorem ConNF.constructMotive_allPermSderiv_forget [Params] {α : Λ} (M : (β : Λ) → β < αMotive β) (H : (β : Λ) → (h : β < α) → Hypothesis (M β h) fun (γ : Λ) (h' : γ < β) => M γ ) {β : Λ} (h : β < α) (ρ : AllPerm α) :
        theorem ConNF.constructMotive_allPermBotSderiv_forget [Params] {α : Λ} (M : (β : Λ) → β < αMotive β) (H : (β : Λ) → (h : β < α) → Hypothesis (M β h) fun (γ : Λ) (h' : γ < β) => M γ ) (ρ : AllPerm α) :
        theorem ConNF.constructMotive_pos_atom_lt_pos [Params] {α : Λ} (M : (β : Λ) → β < αMotive β) (H : (β : Λ) → (h : β < α) → Hypothesis (M β h) fun (γ : Λ) (h' : γ < β) => M γ ) (t : Tangle α) (A : α ) (a : Atom) :
        a (t.support ⇘. A)pos a < pos t
        theorem ConNF.constructMotive_pos_nearLitter_lt_pos [Params] {α : Λ} (M : (β : Λ) → β < αMotive β) (H : (β : Λ) → (h : β < α) → Hypothesis (M β h) fun (γ : Λ) (h' : γ < β) => M γ ) (t : Tangle α) (A : α ) (M✝ : NearLitter) :
        M✝ (t.support ⇘. A)pos M✝ < pos t
        theorem ConNF.constructMotive_smul_fuzz [Params] {α : Λ} (M : (β : Λ) → β < αMotive β) (H : (β : Λ) → (h : β < α) → Hypothesis (M β h) fun (γ : Λ) (h' : γ < β) => M γ ) {β γ : Λ} ( : β < α) ( : γ < α) (hβγ : β γ) (ρ : AllPerm α) (t : Tangle β) :
        theorem ConNF.constructMotive_smul_fuzz_bot [Params] {α : Λ} (M : (β : Λ) → β < αMotive β) (H : (β : Λ) → (h : β < α) → Hypothesis (M β h) fun (γ : Λ) (h' : γ < β) => M γ ) {γ : Λ} ( : γ < α) (ρ : AllPerm α) (t : Tangle ) :
        theorem ConNF.constructMotive_allPerm_of_smul_fuzz [Params] {α : Λ} (M : (β : Λ) → β < αMotive β) (H : (β : Λ) → (h : β < α) → Hypothesis (M β h) fun (γ : Λ) (h' : γ < β) => M γ ) (ρs : {β : Λ} → ( : β < α) → AllPerm β) (π : AllPerm ) :
        (∀ {β γ : Λ} ( : β < α) ( : γ < α) (hδε : β γ) (t : Tangle β), (ρs ) ↘. fuzz hδε t = fuzz hδε (ρs t))(∀ {γ : Λ} ( : γ < α) (t : Tangle ), (ρs ) ↘. fuzz t = fuzz (π t))∃ (ρ : AllPerm α), (∀ (β : Λ) ( : β < α), constructAllPermSderiv M H ρ = ρs ) constructAllPermBotSderiv M H ρ = π
        theorem ConNF.constructMotive_tSet_ext [Params] {α : Λ} (M : (β : Λ) → β < αMotive β) (H : (β : Λ) → (h : β < α) → Hypothesis (M β h) fun (γ : Λ) (h' : γ < β) => M γ ) (β : Λ) ( : β < α) (x y : TSet α) :
        (∀ (z : TSet β), z ∈[] x z ∈[] y)x = y
        theorem ConNF.constructMotive_typedMem_singleton_iff [Params] {α : Λ} (M : (β : Λ) → β < αMotive β) (H : (β : Λ) → (h : β < α) → Hypothesis (M β h) fun (γ : Λ) (h' : γ < β) => M γ ) {β : Λ} ( : β < α) (x y : TSet β) :
        y ∈[] constructSingleton M H x y = x
        def ConNF.constructHypothesis [Params] (α : Λ) (M : (β : Λ) → β < αMotive β) (H : (β : Λ) → (h : β < α) → Hypothesis (M β h) fun (γ : Λ) (h' : γ < β) => M γ ) :
        Equations
        • One or more equations did not get rendered due to their size.
        Instances For