src/HOL/UNITY/PPROD.ML
changeset 10834 a7897aebbffc
parent 10064 1a77667b21ef
child 11220 db536a42dfc5
equal deleted inserted replaced
10833:c0844a30ea4e 10834:a7897aebbffc
   125 \       OK I (%i. lift i (F i)) |]  \
   125 \       OK I (%i. lift i (F i)) |]  \
   126 \    ==> (PLam I F) : X guarantees Y"; 
   126 \    ==> (PLam I F) : X guarantees Y"; 
   127 by (asm_simp_tac (simpset() addsimps [guarantees_JN_I]) 1);
   127 by (asm_simp_tac (simpset() addsimps [guarantees_JN_I]) 1);
   128 qed "guarantees_PLam_I";
   128 qed "guarantees_PLam_I";
   129 
   129 
   130 Goal "Allowed (PLam I F) = (INT i:I. lift i `` Allowed(F i))";
   130 Goal "Allowed (PLam I F) = (INT i:I. lift i ` Allowed(F i))";
   131 by (simp_tac (simpset() addsimps [PLam_def]) 1); 
   131 by (simp_tac (simpset() addsimps [PLam_def]) 1); 
   132 qed "Allowed_PLam";
   132 qed "Allowed_PLam";
   133 Addsimps [Allowed_PLam];
   133 Addsimps [Allowed_PLam];
   134 
   134 
   135 Goal "(PLam I F) : preserves v = (ALL i:I. F i : preserves (v o lift_map i))";
   135 Goal "(PLam I F) : preserves v = (ALL i:I. F i : preserves (v o lift_map i))";