Quot/Examples/SigmaEx.thy
changeset 908 1bf4337919d3
parent 905 51e5cc3793d2
child 912 aa960d16570f
equal deleted inserted replaced
907:e576a97e9a3e 908:1bf4337919d3
   139  (\<forall>l m. hom_e (l, m) = fpar (hom_m m) l m) \<and>
   139  (\<forall>l m. hom_e (l, m) = fpar (hom_m m) l m) \<and>
   140  (\<forall>x a. hom_m (Sig x a) = fsgm (\<lambda>y. hom_o ([(x, y)] \<bullet> a)) (\<lambda>y. [(x, y)] \<bullet> a))
   140  (\<forall>x a. hom_m (Sig x a) = fsgm (\<lambda>y. hom_o ([(x, y)] \<bullet> a)) (\<lambda>y. [(x, y)] \<bullet> a))
   141 )"
   141 )"
   142 apply (lifting tolift)
   142 apply (lifting tolift)
   143 apply (regularize)
   143 apply (regularize)
       
   144 apply (simp)
   144 prefer 2
   145 prefer 2
   145 apply cleaning
   146 apply cleaning
   146 apply simp
   147 apply simp
   147 sorry
   148 sorry
   148 
   149