resolved conflict
authornipkow
Fri, 18 Jan 2019 21:22:46 +0100
changeset 69686 aeceb14f387a
parent 69684 94284d4dab98 (current diff)
parent 69685 32eeb55d4bf3 (diff)
child 69687 b18353d3fe1a
resolved conflict
src/HOL/Analysis/Cartesian_Euclidean_Space.thy
src/HOL/Analysis/Finite_Product_Measure.thy
--- a/src/HOL/Analysis/Cartesian_Euclidean_Space.thy	Thu Jan 17 17:50:01 2019 -0500
+++ b/src/HOL/Analysis/Cartesian_Euclidean_Space.thy	Fri Jan 18 21:22:46 2019 +0100
@@ -2,7 +2,7 @@
    Some material by Jose Divasón, Tim Makarios and L C Paulson
 *)
 
-section%important \<open>Instantiates the finite Cartesian product of Euclidean spaces as a Euclidean space\<close>
+section%important \<open>Finite Cartesian Products of Euclidean Spaces\<close>
 
 theory Cartesian_Euclidean_Space
 imports Cartesian_Space Derivative
--- a/src/HOL/Analysis/Finite_Product_Measure.thy	Thu Jan 17 17:50:01 2019 -0500
+++ b/src/HOL/Analysis/Finite_Product_Measure.thy	Fri Jan 18 21:22:46 2019 +0100
@@ -15,7 +15,7 @@
 lemma case_prod_const: "(\<lambda>(i, j). c) = (\<lambda>_. c)"
   by auto
 
-subsubsection \<open>More about Function restricted by \<^const>\<open>extensional\<close>\<close>
+subsection%unimportant \<open>More about Function restricted by \<^const>\<open>extensional\<close>\<close>
 
 definition
   "merge I J = (\<lambda>(x, y) i. if i \<in> I then x i else if i \<in> J then y i else undefined)"
@@ -111,8 +111,14 @@
 
 subsection \<open>Finite product spaces\<close>
 
+<<<<<<< local
 subsubsection \<open>Products\<close>
 
+||||||| base
+subsubsection%important \<open>Products\<close>
+
+=======
+>>>>>>> other
 definition%important prod_emb where
   "prod_emb I M K X = (\<lambda>x. restrict x K) -` X \<inter> (\<Pi>\<^sub>E i\<in>I. space (M i))"